doc-src/IsarRef/Thy/ZF_Specific.thy
changeset 28761 9ec4482c9201
parent 28760 cbc435f7b16b
child 30168 9a20be5be90b
--- a/doc-src/IsarRef/Thy/ZF_Specific.thy	Thu Nov 13 21:43:46 2008 +0100
+++ b/doc-src/IsarRef/Thy/ZF_Specific.thy	Thu Nov 13 21:45:40 2008 +0100
@@ -16,9 +16,9 @@
   Simplifier setup.
 
   \begin{matharray}{rcl}
-    @{command_def (ZF) "print_tcset"}@{text "\<^sup>*"} & : & \isarkeep{theory~|~proof} \\
-    @{method_def (ZF) typecheck} & : & \isarmeth \\
-    @{attribute_def (ZF) TC} & : & \isaratt \\
+    @{command_def (ZF) "print_tcset"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
+    @{method_def (ZF) typecheck} & : & @{text method} \\
+    @{attribute_def (ZF) TC} & : & @{text attribute} \\
   \end{matharray}
 
   \begin{rail}
@@ -51,10 +51,10 @@
   Coinductive definitions are available in both cases, too.
 
   \begin{matharray}{rcl}
-    @{command_def (ZF) "inductive"} & : & \isartrans{theory}{theory} \\
-    @{command_def (ZF) "coinductive"} & : & \isartrans{theory}{theory} \\
-    @{command_def (ZF) "datatype"} & : & \isartrans{theory}{theory} \\
-    @{command_def (ZF) "codatatype"} & : & \isartrans{theory}{theory} \\
+    @{command_def (ZF) "inductive"} & : & @{text "theory \<rightarrow> theory"} \\
+    @{command_def (ZF) "coinductive"} & : & @{text "theory \<rightarrow> theory"} \\
+    @{command_def (ZF) "datatype"} & : & @{text "theory \<rightarrow> theory"} \\
+    @{command_def (ZF) "codatatype"} & : & @{text "theory \<rightarrow> theory"} \\
   \end{matharray}
 
   \begin{rail}
@@ -104,7 +104,7 @@
 
 text {*
   \begin{matharray}{rcl}
-    @{command_def (ZF) "primrec"} & : & \isartrans{theory}{theory} \\
+    @{command_def (ZF) "primrec"} & : & @{text "theory \<rightarrow> theory"} \\
   \end{matharray}
 
   \begin{rail}
@@ -121,10 +121,10 @@
   ported to Isar.  These should not be used in proper proof texts.
 
   \begin{matharray}{rcl}
-    @{method_def (ZF) case_tac}@{text "\<^sup>*"} & : & \isarmeth \\
-    @{method_def (ZF) induct_tac}@{text "\<^sup>*"} & : & \isarmeth \\
-    @{method_def (ZF) ind_cases}@{text "\<^sup>*"} & : & \isarmeth \\
-    @{command_def (ZF) "inductive_cases"} & : & \isartrans{theory}{theory} \\
+    @{method_def (ZF) case_tac}@{text "\<^sup>*"} & : & @{text method} \\
+    @{method_def (ZF) induct_tac}@{text "\<^sup>*"} & : & @{text method} \\
+    @{method_def (ZF) ind_cases}@{text "\<^sup>*"} & : & @{text method} \\
+    @{command_def (ZF) "inductive_cases"} & : & @{text "theory \<rightarrow> theory"} \\
   \end{matharray}
 
   \begin{rail}