avoid clash of terminology wrt. "semi-automated" in the sense of Isar (e.g. method "rule");
authorwenzelm
Sun, 04 Nov 2012 20:23:26 +0100
changeset 50070 e447ad4d6edd
parent 50069 a10fc2bd3182
child 50071 959548c3b947
avoid clash of terminology wrt. "semi-automated" in the sense of Isar (e.g. method "rule");
src/Doc/IsarRef/Generic.thy
--- a/src/Doc/IsarRef/Generic.thy	Sun Nov 04 20:12:01 2012 +0100
+++ b/src/Doc/IsarRef/Generic.thy	Sun Nov 04 20:23:26 2012 +0100
@@ -1189,7 +1189,7 @@
 *}
 
 
-subsection {* Automated methods *}
+subsection {* Fully automated methods *}
 
 text {*
   \begin{matharray}{rcl}
@@ -1324,7 +1324,7 @@
 *}
 
 
-subsection {* Semi-automated methods *}
+subsection {* Partially automated methods *}
 
 text {* These proof methods may help in situations when the
   fully-automated tools fail.  The result is a simpler subgoal that
@@ -1370,9 +1370,9 @@
     @{index_ML clarify_step_tac: "Proof.context -> int -> tactic"} \\
   \end{matharray}
 
-  These are the primitive tactics behind the (semi)automated proof
-  methods of the Classical Reasoner.  By calling them yourself, you
-  can execute these procedures one step at a time.
+  These are the primitive tactics behind the automated proof methods
+  of the Classical Reasoner.  By calling them yourself, you can
+  execute these procedures one step at a time.
 
   \begin{description}