src/HOL/Bali/DeclConcepts.thy
changeset 23747 b07cff284683
parent 22426 1c38ca2496c4
child 24038 18182c4aec9e
--- a/src/HOL/Bali/DeclConcepts.thy	Wed Jul 11 11:14:51 2007 +0200
+++ b/src/HOL/Bali/DeclConcepts.thy	Wed Jul 11 11:16:34 2007 +0200
@@ -541,7 +541,7 @@
    below
 *)
 
-inductive2
+inductive
   members :: "prog \<Rightarrow> (qtname \<times> memberdecl) \<Rightarrow> qtname \<Rightarrow> bool"
     ("_ \<turnstile> _ member'_of _" [61,61,61] 60)
   for G :: prog
@@ -634,7 +634,7 @@
 
 text {* Static overriding (used during the typecheck of the compiler) *}
 
-inductive2
+inductive
   stat_overridesR :: "prog \<Rightarrow> (qtname \<times> mdecl) \<Rightarrow> (qtname \<times> mdecl) \<Rightarrow> bool"
     ("_ \<turnstile> _ overrides\<^sub>S _" [61,61,61] 60)
   for G :: prog
@@ -653,7 +653,7 @@
 
 text {* Dynamic overriding (used during the typecheck of the compiler) *}
 
-inductive2
+inductive
   overridesR :: "prog \<Rightarrow> (qtname \<times> mdecl) \<Rightarrow> (qtname \<times> mdecl) \<Rightarrow> bool"
     ("_ \<turnstile> _ overrides _" [61,61,61] 60)
   for G :: prog
@@ -784,7 +784,7 @@
 \end{itemize} 
 *} 
 
-inductive2
+inductive
   accessible_fromR :: "prog \<Rightarrow> qtname \<Rightarrow> (qtname \<times> memberdecl) \<Rightarrow> qtname \<Rightarrow> bool"
   and accessible_from :: "prog \<Rightarrow> (qtname \<times> memberdecl) \<Rightarrow> qtname \<Rightarrow> qtname \<Rightarrow> bool"
     ("_ \<turnstile> _ of _ accessible'_from _" [61,61,61,61] 60)
@@ -828,7 +828,7 @@
 "G\<turnstile>Field fn f of C accessible_from accclass"  
  \<rightleftharpoons> "G\<turnstile>(fieldm fn f) of C accessible_from accclass" 
 
-inductive2
+inductive
   dyn_accessible_fromR :: "prog \<Rightarrow> qtname \<Rightarrow> (qtname \<times> memberdecl) \<Rightarrow> qtname \<Rightarrow> bool"
   and dyn_accessible_from' ::  "prog \<Rightarrow> (qtname \<times> memberdecl) \<Rightarrow> qtname \<Rightarrow> qtname \<Rightarrow> bool"
     ("_ \<turnstile> _ in _ dyn'_accessible'_from _" [61,61,61,61] 60)