lsp: changed State_Init notification into a request and removed State_Init_Response;
theory Quickcheck_Nesting_Exampleimports Quickcheck_Nestingbegindatatype x = X "x list"lemma "X a = X b"quickcheck[exhaustive, size = 4, expect = counterexample]oopsend