diff -r 19b47bfac6ef -r 9e7d1c139569 src/Doc/IsarRef/ML_Tactic.thy --- a/src/Doc/IsarRef/ML_Tactic.thy Tue Apr 16 17:54:14 2013 +0200 +++ b/src/Doc/IsarRef/ML_Tactic.thy Thu Apr 18 17:07:01 2013 +0200 @@ -88,12 +88,12 @@ \medskip \begin{tabular}{lll} - @{ML asm_full_simp_tac}~@{text "@{simpset} 1"} & & @{method simp} \\ - @{ML ALLGOALS}~(@{ML asm_full_simp_tac}~@{text "@{simpset}"}) & & @{method simp_all} \\[0.5ex] - @{ML simp_tac}~@{text "@{simpset} 1"} & & @{method simp}~@{text "(no_asm)"} \\ - @{ML asm_simp_tac}~@{text "@{simpset} 1"} & & @{method simp}~@{text "(no_asm_simp)"} \\ - @{ML full_simp_tac}~@{text "@{simpset} 1"} & & @{method simp}~@{text "(no_asm_use)"} \\ - @{ML asm_lr_simp_tac}~@{text "@{simpset} 1"} & & @{method simp}~@{text "(asm_lr)"} \\ + @{ML asm_full_simp_tac}~@{text "@{context} 1"} & & @{method simp} \\ + @{ML ALLGOALS}~(@{ML asm_full_simp_tac}~@{text "@{context}"}) & & @{method simp_all} \\[0.5ex] + @{ML simp_tac}~@{text "@{context} 1"} & & @{method simp}~@{text "(no_asm)"} \\ + @{ML asm_simp_tac}~@{text "@{context} 1"} & & @{method simp}~@{text "(no_asm_simp)"} \\ + @{ML full_simp_tac}~@{text "@{context} 1"} & & @{method simp}~@{text "(no_asm_use)"} \\ + @{ML asm_lr_simp_tac}~@{text "@{context} 1"} & & @{method simp}~@{text "(asm_lr)"} \\ \end{tabular} \medskip *}