src/HOL/IMP/Live_True.thy
changeset 68484 59793df7f853
parent 67406 23307fd33906
child 68776 403dd13cf6e9
--- a/src/HOL/IMP/Live_True.thy	Fri Jun 22 18:31:50 2018 +0200
+++ b/src/HOL/IMP/Live_True.thy	Fri Jun 22 20:31:49 2018 +0200
@@ -115,7 +115,7 @@
 qed auto
 
 text\<open>Make @{const L} executable by replacing @{const lfp} with the @{const
-while} combinator from theory @{theory While_Combinator}. The @{const while}
+while} combinator from theory @{theory "HOL-Library.While_Combinator"}. The @{const while}
 combinator obeys the recursion equation
 @{thm[display] While_Combinator.while_unfold[no_vars]}
 and is thus executable.\<close>