(* Title: HOL/Induct/Com.thy Author: Lawrence C Paulson, Cambridge University Computer Laboratory Copyright 1997 University of Cambridge Example of Mutual Induction via Iteratived Inductive Definitions: Commands *) section‹Mutual Induction via Iteratived Inductive Definitions› theory Com imports Main begin typedecl loc type_synonym state = "loc => nat"